aboutsummaryrefslogtreecommitdiffstats
path: root/src/Verilog/VerilogAST.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Verilog/VerilogAST.v')
-rw-r--r--src/Verilog/VerilogAST.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/Verilog/VerilogAST.v b/src/Verilog/VerilogAST.v
index 5886652..8bb8ba8 100644
--- a/src/Verilog/VerilogAST.v
+++ b/src/Verilog/VerilogAST.v
@@ -22,7 +22,8 @@ Structures.OrderedTypeEx
FSets.FMapList
Program.Basics
PeanoNat.
-From CoqUp.Common Require Import Helper Tactics Show.
+
+From coqup.common Require Import Helper Tactics Show.
Import ListNotations.
@@ -32,8 +33,7 @@ Inductive value : Type :=
| VBool (b : bool)
| VArray (l : list value).
-Inductive literal : Type :=
-| LitArray (l : list bool).
+Inductive literal : Type := LitArray (l : list bool).
Definition cons_value (a b : value) : value :=
match a, b with