tuned
authorhaftmann
Mon, 01 Jun 2015 18:59:19 +0200
changeset 60337 c7ca6bb006b0
parent 60336 f0b2457bf68e
child 60338 a808b57d5b0d
tuned
src/Pure/Isar/class.ML
src/Pure/Isar/generic_target.ML
--- a/src/Pure/Isar/class.ML	Mon Jun 01 18:07:36 2015 +0200
+++ b/src/Pure/Isar/class.ML	Mon Jun 01 18:59:19 2015 +0200
@@ -336,7 +336,7 @@
     val rhs2 = Morphism.term phi2 rhs;
   in n1 = n2 andalso Term.aconv_untyped (rhs1, rhs2) end;
 
-fun target_const class phi0 prmode ((b, _), rhs) =
+fun target_const class phi0 prmode (b, rhs) =
   let
     val guess_identity = guess_morphism_identity (b, rhs) Morphism.identity;
     val guess_canonical = guess_morphism_identity (b, rhs) phi0;
@@ -404,7 +404,7 @@
     val dangling_params = map (Morphism.term phi) (uncurry append (dangling_params_for lthy class params));
   in
     lthy
-    |> target_const class phi Syntax.mode_default ((b, mx), lhs)
+    |> target_const class phi Syntax.mode_default (b, lhs)
     |> Local_Theory.raw_theory (canonical_const class phi dangling_params
          ((Morphism.binding phi b, if null dangling_params then mx else NoSyn), Morphism.term phi lhs))
     |> Generic_Target.standard_const (fn (this, other) => other <> 0 andalso this <> other)
@@ -418,7 +418,7 @@
     val dangling_term_params = map (Morphism.term phi) (snd (dangling_params_for lthy class params));
   in
     lthy
-    |> target_const class phi prmode ((b, mx), lhs)
+    |> target_const class phi prmode (b, lhs)
     |> Local_Theory.raw_theory (canonical_abbrev class phi prmode dangling_term_params
          ((Morphism.binding phi b, if null dangling_term_params then mx else NoSyn), rhs'))
     |> Generic_Target.standard_const (fn (this, other) => other <> 0 andalso this <> other)
--- a/src/Pure/Isar/generic_target.ML	Mon Jun 01 18:07:36 2015 +0200
+++ b/src/Pure/Isar/generic_target.ML	Mon Jun 01 18:59:19 2015 +0200
@@ -27,9 +27,9 @@
       (Attrib.binding * (thm list * Token.src list) list) list -> local_theory -> local_theory) ->
     string -> (Attrib.binding * (thm list * Token.src list) list) list -> local_theory ->
     (string * thm list) list * local_theory
-  val abbrev: (string * bool -> binding * mixfix -> term ->
+  val abbrev: (Syntax.mode -> binding * mixfix -> term ->
       term list * term list -> local_theory -> local_theory) ->
-    string * bool -> (binding * mixfix) * term -> local_theory -> (term * term) * local_theory
+    Syntax.mode -> (binding * mixfix) * term -> local_theory -> (term * term) * local_theory
 
   (*theory operations*)
   val theory_foundation: ((binding * typ) * mixfix) * (binding * term) ->