src/HOL/Mutabelle/Mutabelle.thy
changeset 38864 4abe644fcea5
parent 38795 848be46708dc
child 39557 fe5722fce758
--- a/src/HOL/Mutabelle/Mutabelle.thy	Sat Aug 28 20:24:40 2010 +0800
+++ b/src/HOL/Mutabelle/Mutabelle.thy	Sat Aug 28 16:14:32 2010 +0200
@@ -4,7 +4,7 @@
 begin
 
 ML {*
-val comms = [@{const_name "op ="}, @{const_name HOL.disj}, @{const_name HOL.conj}];
+val comms = [@{const_name HOL.eq}, @{const_name HOL.disj}, @{const_name HOL.conj}];
 
 val forbidden =
  [(@{const_name Power.power}, "'a"),