aboutsummaryrefslogtreecommitdiffstats
path: root/src/Extraction/Extraction.v
blob: c4248cb7e5e43e572c390192698d83bce713ea0e (plain)
1
2
3
4
5
6
7
8
Require CoqUp.Verilog.VerilogAST.

Require Import ExtrOcamlBasic.
Require Import ExtrOcamlString.

Cd "src/Extraction".
Separate Extraction
         VerilogAST.nat_to_value VerilogAST.value_to_nat VerilogAST.verilog VerilogAST.verilog_example.