new datatype is too slow on the huge datatypes (at least the mutual ones) -- use 'old_datatype' instead
authorblanchet
Fri, 12 Sep 2014 17:30:05 +0200
changeset 58330 a016c42d136d
parent 58329 a31404ec7414
child 58331 054e9a9fccad
new datatype is too slow on the huge datatypes (at least the mutual ones) -- use 'old_datatype' instead
src/HOL/Datatype_Examples/Brackin.thy
src/HOL/Datatype_Examples/Instructions.thy
src/HOL/Datatype_Examples/SML.thy
src/HOL/Datatype_Examples/Verilog.thy
--- a/src/HOL/Datatype_Examples/Brackin.thy	Fri Sep 12 16:42:36 2014 +0200
+++ b/src/HOL/Datatype_Examples/Brackin.thy	Fri Sep 12 17:30:05 2014 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Datatype_Benchmark/Brackin.thy
+(*  Title:      HOL/Datatype_Examples/Brackin.thy
 
 A couple of datatypes from Steve Brackin's work.
 *)
--- a/src/HOL/Datatype_Examples/Instructions.thy	Fri Sep 12 16:42:36 2014 +0200
+++ b/src/HOL/Datatype_Examples/Instructions.thy	Fri Sep 12 17:30:05 2014 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Datatype_Benchmark/Instructions.thy
+(*  Title:      HOL/Datatype_Examples/Instructions.thy
 
 Example from Konrad: 68000 instruction set.
 *)
@@ -59,7 +59,7 @@
 | pcdisp nat
 | pcindex nat DataOrAddressRegister Size
 
-datatype M68kInstruction =
+old_datatype M68kInstruction =
   ABCD AddressingMode AddressingMode
 | ADD Size AddressingMode AddressingMode
 | ADDA Size AddressingMode AddressRegister
--- a/src/HOL/Datatype_Examples/SML.thy	Fri Sep 12 16:42:36 2014 +0200
+++ b/src/HOL/Datatype_Examples/SML.thy	Fri Sep 12 17:30:05 2014 +0200
@@ -1,4 +1,4 @@
-(*  Title:      HOL/Datatype_Benchmark/SML.thy
+(*  Title:      HOL/Datatype_Examples/SML.thy
 
 Example from Myra: part of the syntax of SML.
 *)
@@ -32,7 +32,7 @@
 datatype
   'a long = BASE 'a | QUALIFIED strid "'a long"
 
-datatype
+old_datatype
    atpat_e = WILDCARDatpat_e
            | SCONatpat_e scon
            | VARatpat_e var
--- a/src/HOL/Datatype_Examples/Verilog.thy	Fri Sep 12 16:42:36 2014 +0200
+++ b/src/HOL/Datatype_Examples/Verilog.thy	Fri Sep 12 17:30:05 2014 +0200
@@ -1,11 +1,11 @@
-(*  Title:      HOL/Datatype_Benchmark/Verilog.thy
+(*  Title:      HOL/Datatype_Examples/Verilog.thy
 
 Example from Daryl: a Verilog grammar.
 *)
 
 theory Verilog imports Main begin
 
-datatype
+old_datatype
   Source_text
      = module string "string list" "Module_item list"
      | Source_textMeta string