Quot/quotient_term.ML
author Cezary Kaliszyk <kaliszyk@in.tum.de>
Wed, 13 Jan 2010 16:23:32 +0100
changeset 865 5c6d76c3ba5c
parent 858 bb012513fb39
child 867 9e247b9505f0
permissions -rw-r--r--
Put relation_error as a separate function.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     1
signature QUOTIENT_TERM =
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
     2
sig
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
     3
  exception LIFT_MATCH of string
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
     4
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
     5
  datatype flag = absF | repF
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
     6
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
     7
  val absrep_fun: flag -> Proof.context -> typ * typ -> term
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
     8
  val absrep_fun_chk: flag -> Proof.context -> typ * typ -> term
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
     9
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    10
  val equiv_relation: Proof.context -> typ * typ -> term
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    11
  val equiv_relation_chk: Proof.context -> typ * typ -> term
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
    12
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    13
  val regularize_trm: Proof.context -> term * term -> term
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    14
  val regularize_trm_chk: Proof.context -> term * term -> term
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    15
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    16
  val inj_repabs_trm: Proof.context -> term * term -> term
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    17
  val inj_repabs_trm_chk: Proof.context -> term * term -> term
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    18
end;
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    19
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    20
structure Quotient_Term: QUOTIENT_TERM =
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    21
struct
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
    22
762
baac4639ecef avoided global "open"s - replaced by local "open"s
Christian Urban <urbanc@in.tum.de>
parents: 761
diff changeset
    23
open Quotient_Info;
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    24
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    25
exception LIFT_MATCH of string
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    26
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
    27
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
    28
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
    29
(*** Aggregate Rep/Abs Function ***)
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
    30
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
    31
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    32
(* The flag repF is for types in negative position; absF is for types 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    33
   in positive position. Because of this, function types need to be   
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    34
   treated specially, since there the polarity changes.               
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    35
*)
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    36
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    37
datatype flag = absF | repF
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    38
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    39
fun negF absF = repF
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    40
  | negF repF = absF
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    41
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    42
fun is_identity (Const (@{const_name "id"}, _)) = true
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    43
  | is_identity _ = false
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    44
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    45
fun mk_identity ty = Const (@{const_name "id"}, ty --> ty)
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    46
807
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
    47
fun mk_fun_compose flag (trm1, trm2) = 
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    48
  case flag of
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    49
    absF => Const (@{const_name "comp"}, dummyT) $ trm1 $ trm2
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    50
  | repF => Const (@{const_name "comp"}, dummyT) $ trm2 $ trm1
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    51
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    52
fun get_mapfun ctxt s =
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    53
let
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
    54
  val thy = ProofContext.theory_of ctxt
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    55
  val exc = LIFT_MATCH ("No map function for type " ^ quote s ^ " found.")
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    56
  val mapfun = #mapfun (maps_lookup thy s) handle NotFound => raise exc
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    57
in
784
da75568e7f12 renamed some fields in the info records
Christian Urban <urbanc@in.tum.de>
parents: 783
diff changeset
    58
  Const (mapfun, dummyT)
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    59
end
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    60
800
71225f4a4635 some slight tuning
Christian Urban <urbanc@in.tum.de>
parents: 797
diff changeset
    61
(* makes a Free out of a TVar *)
71225f4a4635 some slight tuning
Christian Urban <urbanc@in.tum.de>
parents: 797
diff changeset
    62
fun mk_Free (TVar ((x, i), _)) = Free (unprefix "'" x ^ string_of_int i, dummyT)
71225f4a4635 some slight tuning
Christian Urban <urbanc@in.tum.de>
parents: 797
diff changeset
    63
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    64
(* produces an aggregate map function for the       
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    65
   rty-part of a quotient definition; abstracts     
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    66
   over all variables listed in vs (these variables 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    67
   correspond to the type variables in rty)         
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    68
                                                    
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    69
   for example for: (?'a list * ?'b)                
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    70
   it produces:     %a b. prod_map (map a) b 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    71
*)
803
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
    72
fun mk_mapfun ctxt vs rty =
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    73
let
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    74
  val vs' = map (mk_Free) vs
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    75
803
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
    76
  fun mk_mapfun_aux rty =
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
    77
    case rty of
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
    78
      TVar _ => mk_Free rty
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
    79
    | Type (_, []) => mk_identity rty
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    80
    | Type (s, tys) => list_comb (get_mapfun ctxt s, map mk_mapfun_aux tys)
804
Christian Urban <urbanc@in.tum.de>
parents: 803
diff changeset
    81
    | _ => raise LIFT_MATCH ("mk_mapfun (default)")
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    82
in
803
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
    83
  fold_rev Term.lambda vs' (mk_mapfun_aux rty)
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    84
end
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    85
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    86
(* looks up the (varified) rty and qty for 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    87
   a quotient definition                   
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    88
*)
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    89
fun get_rty_qty ctxt s =
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
    90
let
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
    91
  val thy = ProofContext.theory_of ctxt
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
    92
  val exc = LIFT_MATCH ("No quotient type " ^ quote s ^ " found.")
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    93
  val qdata = (quotdata_lookup thy s) handle NotFound => raise exc
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    94
in
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    95
  (#rtyp qdata, #qtyp qdata)
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    96
end
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
    97
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    98
(* takes two type-environments and looks    
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
    99
   up in both of them the variable v, which 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   100
   must be listed in the environment        
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   101
*)
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   102
fun double_lookup rtyenv qtyenv v =
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   103
let
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   104
  val v' = fst (dest_TVar v)
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   105
in
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   106
  (snd (the (Vartab.lookup rtyenv v')), snd (the (Vartab.lookup qtyenv v')))
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   107
end
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   108
832
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   109
(* matches a type pattern with a type *)
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   110
fun match ctxt err ty_pat ty =
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   111
let
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   112
  val thy = ProofContext.theory_of ctxt
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   113
in
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   114
  Sign.typ_match thy (ty_pat, ty) Vartab.empty
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   115
  handle MATCH_TYPE => err ctxt ty_pat ty
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   116
end
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   117
800
71225f4a4635 some slight tuning
Christian Urban <urbanc@in.tum.de>
parents: 797
diff changeset
   118
(* produces the rep or abs constant for a qty *)
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   119
fun absrep_const flag ctxt qty_str =
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   120
let
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   121
  val thy = ProofContext.theory_of ctxt
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   122
  val qty_name = Long_Name.base_name qty_str
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   123
in
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   124
  case flag of
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   125
    absF => Const (Sign.full_bname thy ("abs_" ^ qty_name), dummyT)
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   126
  | repF => Const (Sign.full_bname thy ("rep_" ^ qty_name), dummyT)
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   127
end
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   128
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   129
fun absrep_match_err ctxt ty_pat ty =
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   130
let
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   131
  val ty_pat_str = Syntax.string_of_typ ctxt ty_pat
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   132
  val ty_str = Syntax.string_of_typ ctxt ty 
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   133
in
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   134
  raise LIFT_MATCH (space_implode " " 
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   135
    ["absrep_fun (Types ", quote ty_pat_str, "and", quote ty_str, " do not match.)"])
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   136
end
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   137
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   138
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   139
(** generation of an aggregate absrep function **)
791
fb4bfbb1a291 commeted the absrep function
Christian Urban <urbanc@in.tum.de>
parents: 790
diff changeset
   140
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   141
(* - In case of equal types we just return the identity.           
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   142
     
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   143
   - In case of TFrees we also return the identity.
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   144
                                                             
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   145
   - In case of function types we recurse taking   
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   146
     the polarity change into account.              
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   147
                                                                   
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   148
   - If the type constructors are equal, we recurse for the        
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   149
     arguments and build the appropriate map function.             
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   150
                                                                   
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   151
   - If the type constructors are unequal, there must be an        
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   152
     instance of quotient types:         
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   153
                          
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   154
       - we first look up the corresponding rty_pat and qty_pat    
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   155
         from the quotient definition; the arguments of qty_pat    
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   156
         must be some distinct TVars                               
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   157
       - we then match the rty_pat with rty and qty_pat with qty;  
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   158
         if matching fails the types do not correspond -> error                  
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   159
       - the matching produces two environments; we look up the    
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   160
         assignments for the qty_pat variables and recurse on the  
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   161
         assignments                                               
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   162
       - we prefix the aggregate map function for the rty_pat,     
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   163
         which is an abstraction over all type variables           
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   164
       - finally we compose the result with the appropriate        
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   165
         absrep function in case at least one argument produced
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   166
         a non-identity function /
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   167
         otherwise we just return the appropriate absrep
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   168
         function                                          
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   169
                                                                   
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   170
     The composition is necessary for types like                   
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   171
                                                                 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   172
        ('a list) list / ('a foo) foo                              
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   173
                                                                 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   174
     The matching is necessary for types like                      
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   175
                                                                 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   176
        ('a * 'a) list / 'a bar   
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   177
858
Christian Urban <urbanc@in.tum.de>
parents: 856
diff changeset
   178
     The test is necessary in order to eliminate superfluous
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   179
     identity maps.                                 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   180
*)  
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   181
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   182
fun absrep_fun flag ctxt (rty, qty) =
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   183
  if rty = qty  
803
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
   184
  then mk_identity rty
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   185
  else
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   186
    case (rty, qty) of
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   187
      (Type ("fun", [ty1, ty2]), Type ("fun", [ty1', ty2'])) =>
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   188
        let
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   189
          val arg1 = absrep_fun (negF flag) ctxt (ty1, ty1')
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   190
          val arg2 = absrep_fun flag ctxt (ty2, ty2')
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   191
        in
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   192
          list_comb (get_mapfun ctxt "fun", [arg1, arg2])
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   193
        end
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   194
    | (Type (s, tys), Type (s', tys')) =>
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   195
        if s = s'
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   196
        then 
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   197
           let
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   198
             val args = map (absrep_fun flag ctxt) (tys ~~ tys')
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   199
           in
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   200
             list_comb (get_mapfun ctxt s, args)
832
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   201
           end 
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   202
        else
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   203
           let
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   204
             val (rty_pat, qty_pat as Type (_, vs)) = get_rty_qty ctxt s'
832
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   205
             val rtyenv = match ctxt absrep_match_err rty_pat rty
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   206
             val qtyenv = match ctxt absrep_match_err qty_pat qty
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   207
             val args_aux = map (double_lookup rtyenv qtyenv) vs
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   208
             val args = map (absrep_fun flag ctxt) args_aux
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   209
             val map_fun = mk_mapfun ctxt vs rty_pat       
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   210
             val result = list_comb (map_fun, args) 
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   211
           in
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   212
             if forall is_identity args
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   213
             then absrep_const flag ctxt s'
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   214
             else mk_fun_compose flag (absrep_const flag ctxt s', result)
830
89d772dae4d4 New_relations, all works again including concat examples.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 826
diff changeset
   215
           end
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   216
    | (TFree x, TFree x') =>
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   217
        if x = x'
803
6f6ee78c7357 a slight change to abs/rep generation
Christian Urban <urbanc@in.tum.de>
parents: 801
diff changeset
   218
        then mk_identity rty
790
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   219
        else raise (LIFT_MATCH "absrep_fun (frees)")
3a48ffcf0f9a generalised absrep function; needs consolidation
Christian Urban <urbanc@in.tum.de>
parents: 786
diff changeset
   220
    | (TVar _, TVar _) => raise (LIFT_MATCH "absrep_fun (vars)")
791
fb4bfbb1a291 commeted the absrep function
Christian Urban <urbanc@in.tum.de>
parents: 790
diff changeset
   221
    | _ => raise (LIFT_MATCH "absrep_fun (default)")
774
b4ffb8826105 moved get_fun into quotient_term; this simplifies the overall including structure of the package
Christian Urban <urbanc@in.tum.de>
parents: 762
diff changeset
   222
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   223
fun absrep_fun_chk flag ctxt (rty, qty) =
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   224
  absrep_fun flag ctxt (rty, qty)
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   225
  |> Syntax.check_term ctxt
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   226
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   227
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   228
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   229
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   230
(*** Aggregate Equivalence Relation ***)
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   231
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   232
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   233
(* works very similar to the absrep generation,
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   234
   except there is no need for polarities
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   235
*)
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   236
783
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   237
(* instantiates TVars so that the term is of type ty *)
792
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   238
fun force_typ ctxt trm ty =
783
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   239
let
792
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   240
  val thy = ProofContext.theory_of ctxt 
783
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   241
  val trm_ty = fastype_of trm
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   242
  val ty_inst = Sign.typ_match thy (trm_ty, ty) Vartab.empty
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   243
in
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   244
  map_types (Envir.subst_type ty_inst) trm
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   245
end
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   246
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   247
fun is_eq (Const (@{const_name "op ="}, _)) = true
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   248
  | is_eq _ = false
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   249
825
970e86082cd7 Modifictaions for new_relation.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 808
diff changeset
   250
fun mk_rel_compose (trm1, trm2) =
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   251
  Const (@{const_name "rel_conj"}, dummyT) $ trm1 $ trm2
807
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   252
792
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   253
fun get_relmap ctxt s =
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   254
let
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   255
  val thy = ProofContext.theory_of ctxt
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   256
  val exc =  LIFT_MATCH ("get_relmap (no relation map function found for type " ^ s ^ ")") 
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   257
  val relmap =  #relmap (maps_lookup thy s) handle NotFound => raise exc
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   258
in
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   259
  Const (relmap, dummyT)
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   260
end
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   261
807
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   262
fun mk_relmap ctxt vs rty =
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   263
let
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   264
  val vs' = map (mk_Free) vs
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   265
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   266
  fun mk_relmap_aux rty =
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   267
    case rty of
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   268
      TVar _ => mk_Free rty
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   269
    | Type (_, []) => HOLogic.eq_const rty
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   270
    | Type (s, tys) => list_comb (get_relmap ctxt s, map mk_relmap_aux tys)
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   271
    | _ => raise LIFT_MATCH ("mk_relmap (default)")
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   272
in
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   273
  fold_rev Term.lambda vs' (mk_relmap_aux rty)
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   274
end
a5495a323b49 added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest)
Christian Urban <urbanc@in.tum.de>
parents: 804
diff changeset
   275
792
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   276
fun get_equiv_rel ctxt s =
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   277
let
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   278
  val thy = ProofContext.theory_of ctxt
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   279
  val exc = LIFT_MATCH ("get_quotdata (no quotient found for type " ^ s ^ ")") 
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   280
in
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   281
  #equiv_rel (quotdata_lookup thy s) handle NotFound => raise exc
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   282
end
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   283
808
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   284
fun equiv_match_err ctxt ty_pat ty =
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   285
let
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   286
  val ty_pat_str = Syntax.string_of_typ ctxt ty_pat
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   287
  val ty_str = Syntax.string_of_typ ctxt ty 
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   288
in
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   289
  raise LIFT_MATCH (space_implode " " 
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   290
    ["equiv_relation (Types ", quote ty_pat_str, "and", quote ty_str, " do not match.)"])
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   291
end
90bde96f5dd1 proper handling of error messages (code copy - maybe this can be avoided)
Christian Urban <urbanc@in.tum.de>
parents: 807
diff changeset
   292
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   293
(* builds the aggregate equivalence relation 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   294
   that will be the argument of Respects     
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   295
*)
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   296
fun equiv_relation ctxt (rty, qty) =
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   297
  if rty = qty
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   298
  then HOLogic.eq_const rty
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   299
  else
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   300
    case (rty, qty) of
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   301
      (Type (s, tys), Type (s', tys')) =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   302
       if s = s' 
761
e2ac18492c68 small tuning
Christian Urban <urbanc@in.tum.de>
parents: 760
diff changeset
   303
       then 
e2ac18492c68 small tuning
Christian Urban <urbanc@in.tum.de>
parents: 760
diff changeset
   304
         let
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   305
           val args = map (equiv_relation ctxt) (tys ~~ tys')
761
e2ac18492c68 small tuning
Christian Urban <urbanc@in.tum.de>
parents: 760
diff changeset
   306
         in
792
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   307
           list_comb (get_relmap ctxt s, args) 
761
e2ac18492c68 small tuning
Christian Urban <urbanc@in.tum.de>
parents: 760
diff changeset
   308
         end  
e2ac18492c68 small tuning
Christian Urban <urbanc@in.tum.de>
parents: 760
diff changeset
   309
       else 
784
da75568e7f12 renamed some fields in the info records
Christian Urban <urbanc@in.tum.de>
parents: 783
diff changeset
   310
         let
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   311
           val (rty_pat, qty_pat as Type (_, vs)) = get_rty_qty ctxt s'
832
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   312
           val rtyenv = match ctxt equiv_match_err rty_pat rty
b3bb2bad952f introduced separate match function
Christian Urban <urbanc@in.tum.de>
parents: 831
diff changeset
   313
           val qtyenv = match ctxt equiv_match_err qty_pat qty
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   314
           val args_aux = map (double_lookup rtyenv qtyenv) vs 
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   315
           val args = map (equiv_relation ctxt) args_aux
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   316
           val rel_map = mk_relmap ctxt vs rty_pat       
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   317
           val result = list_comb (rel_map, args)
792
Christian Urban <urbanc@in.tum.de>
parents: 791
diff changeset
   318
           val eqv_rel = get_equiv_rel ctxt s'
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   319
           val eqv_rel' = force_typ ctxt eqv_rel ([rty, rty] ---> @{typ bool})
761
e2ac18492c68 small tuning
Christian Urban <urbanc@in.tum.de>
parents: 760
diff changeset
   320
         in
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   321
           if forall is_eq args 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   322
           then eqv_rel'
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   323
           else mk_rel_compose (result, eqv_rel')
761
e2ac18492c68 small tuning
Christian Urban <urbanc@in.tum.de>
parents: 760
diff changeset
   324
         end
783
06e17083e90b modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants
Christian Urban <urbanc@in.tum.de>
parents: 782
diff changeset
   325
      | _ => HOLogic.eq_const rty
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   326
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   327
fun equiv_relation_chk ctxt (rty, qty) =
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   328
  equiv_relation ctxt (rty, qty)
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   329
  |> Syntax.check_term ctxt
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   330
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   331
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   332
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   333
(*** Regularization ***)
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   334
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   335
(* Regularizing an rtrm means:
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   336
 
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   337
 - Quantifiers over types that need lifting are replaced 
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   338
   by bounded quantifiers, for example:
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   339
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   340
      All P  ----> All (Respects R) P
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   341
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   342
   where the aggregate relation R is given by the rty and qty;
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   343
 
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   344
 - Abstractions over types that need lifting are replaced
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   345
   by bounded abstractions, for example:
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   346
      
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   347
      %x. P  ----> Ball (Respects R) %x. P
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   348
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   349
 - Equalities over types that need lifting are replaced by
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   350
   corresponding equivalence relations, for example:
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   351
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   352
      A = B  ----> R A B
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   353
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
   354
   or
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   355
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   356
      A = B  ----> (R ===> R) A B
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
   357
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   358
   for more complicated types of A and B
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   359
*)
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   360
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   361
val mk_babs = Const (@{const_name Babs}, dummyT)
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   362
val mk_ball = Const (@{const_name Ball}, dummyT)
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   363
val mk_bex  = Const (@{const_name Bex}, dummyT)
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   364
val mk_resp = Const (@{const_name Respects}, dummyT)
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   365
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   366
(* - applies f to the subterm of an abstraction, 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   367
     otherwise to the given term,                
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   368
   - used by regularize, therefore abstracted    
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   369
     variables do not have to be treated specially 
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   370
*)
775
Christian Urban <urbanc@in.tum.de>
parents: 774
diff changeset
   371
fun apply_subt f (trm1, trm2) =
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   372
  case (trm1, trm2) of
775
Christian Urban <urbanc@in.tum.de>
parents: 774
diff changeset
   373
    (Abs (x, T, t), Abs (_ , _, t')) => Abs (x, T, f (t, t'))
Christian Urban <urbanc@in.tum.de>
parents: 774
diff changeset
   374
  | _ => f (trm1, trm2)
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   375
865
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   376
fun relation_error ctxt r1 r2 =
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   377
let
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   378
  val r1s = Syntax.string_of_term ctxt r1
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   379
  val r2s = Syntax.string_of_term ctxt r2
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   380
  val r1t = Syntax.string_of_typ ctxt (fastype_of r1)
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   381
  val r2t = Syntax.string_of_typ ctxt (fastype_of r2)
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   382
in
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   383
  raise LIFT_MATCH ("regularise (relation mismatch)\n[" ^
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   384
  r1s ^ " :: " ^ r1t ^ "]\n[" ^ r2s ^ " :: " ^ r2t ^ "]")
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   385
end
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   386
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   387
(* the major type of All and Ex quantifiers *)
853
3fd1365f5729 More indenting, bracket removing and comment restructuring.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 849
diff changeset
   388
fun qnt_typ ty = domain_type (domain_type ty)
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   389
856
Christian Urban <urbanc@in.tum.de>
parents: 854 853
diff changeset
   390
(* produces a regularized version of rtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   391
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   392
   - the result might contain dummyTs           
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   393
854
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   394
   - for regularisation we do not need any      
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   395
     special treatment of bound variables       
5961edda27d7 absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 836
diff changeset
   396
*)
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   397
fun regularize_trm ctxt (rtrm, qtrm) =
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   398
  case (rtrm, qtrm) of
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   399
    (Abs (x, ty, t), Abs (_, ty', t')) =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   400
       let
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   401
         val subtrm = Abs(x, ty, regularize_trm ctxt (t, t'))
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   402
       in
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   403
         if ty = ty' then subtrm
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   404
         else mk_babs $ (mk_resp $ equiv_relation ctxt (ty, ty')) $ subtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   405
       end
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   406
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   407
  | (Const (@{const_name "All"}, ty) $ t, Const (@{const_name "All"}, ty') $ t') =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   408
       let
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   409
         val subtrm = apply_subt (regularize_trm ctxt) (t, t')
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   410
       in
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   411
         if ty = ty' then Const (@{const_name "All"}, ty) $ subtrm
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   412
         else mk_ball $ (mk_resp $ equiv_relation ctxt (qnt_typ ty, qnt_typ ty')) $ subtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   413
       end
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   414
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   415
  | (Const (@{const_name "Ex"}, ty) $ t, Const (@{const_name "Ex"}, ty') $ t') =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   416
       let
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   417
         val subtrm = apply_subt (regularize_trm ctxt) (t, t')
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   418
       in
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   419
         if ty = ty' then Const (@{const_name "Ex"}, ty) $ subtrm
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   420
         else mk_bex $ (mk_resp $ equiv_relation ctxt (qnt_typ ty, qnt_typ ty')) $ subtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   421
       end
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   422
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   423
  | (* equalities need to be replaced by appropriate equivalence relations *) 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   424
    (Const (@{const_name "op ="}, ty), Const (@{const_name "op ="}, ty')) =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   425
         if ty = ty' then rtrm
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   426
         else equiv_relation ctxt (domain_type ty, domain_type ty') 
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   427
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   428
  | (* in this case we just check whether the given equivalence relation is correct *) 
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   429
    (rel, Const (@{const_name "op ="}, ty')) =>
865
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   430
       let
785
Christian Urban <urbanc@in.tum.de>
parents: 784
diff changeset
   431
         val rel_ty = fastype_of rel
831
224909b9399f removed obsolete equiv_relation and rnamed new_equiv_relation
Christian Urban <urbanc@in.tum.de>
parents: 830
diff changeset
   432
         val rel' = equiv_relation_chk ctxt (domain_type rel_ty, domain_type ty') 
865
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   433
       in
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   434
         if rel' aconv rel then rtrm else relation_error ctxt rel rel'
5c6d76c3ba5c Put relation_error as a separate function.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 858
diff changeset
   435
       end
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   436
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   437
  | (_, Const _) =>
835
c4fa87dd0208 Fix for testing matching constants in regularize.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 834
diff changeset
   438
       let
c4fa87dd0208 Fix for testing matching constants in regularize.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 834
diff changeset
   439
         val thy = ProofContext.theory_of ctxt
836
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   440
         fun matches_typ T T' =
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   441
           case (T, T') of
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   442
             (TFree _, TFree _) => true
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   443
           | (TVar _, TVar _) => true
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   444
           | (Type (s, tys), Type (s', tys')) => (
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   445
               (s = s' andalso tys = tys') orelse
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   446
               (* 'andalso' is buildin syntax so it needs to be expanded *)
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   447
               (fold (fn x => fn y => x andalso y) (map2 matches_typ tys tys') (s = s')
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   448
                handle UnequalLengths => false
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   449
               ) orelse
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   450
               let
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   451
                 val rty = #rtyp (Quotient_Info.quotdata_lookup thy s')
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   452
               in
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   453
                 Sign.typ_instance thy (T, rty)
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   454
               end
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   455
               handle Not_found => false (* raised by quotdata_lookup *)
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   456
             )
c2501b2b262a removed quotdata_lookup_type
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 835
diff changeset
   457
           | _ => false
835
c4fa87dd0208 Fix for testing matching constants in regularize.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 834
diff changeset
   458
         fun same_const (Const (s, T)) (Const (s', T')) = (s = s') andalso matches_typ T T'
c4fa87dd0208 Fix for testing matching constants in regularize.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 834
diff changeset
   459
           | same_const _ _ = false
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   460
       in
835
c4fa87dd0208 Fix for testing matching constants in regularize.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 834
diff changeset
   461
         if same_const rtrm qtrm then rtrm
c4fa87dd0208 Fix for testing matching constants in regularize.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 834
diff changeset
   462
         else
c4fa87dd0208 Fix for testing matching constants in regularize.
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 834
diff changeset
   463
           let
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   464
             val qtrm_str = Syntax.string_of_term ctxt qtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   465
             val exc1 = LIFT_MATCH ("regularize (constant " ^ qtrm_str ^ " not found)")
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   466
             val exc2 = LIFT_MATCH ("regularize (constant " ^ qtrm_str ^ " mismatch)")
785
Christian Urban <urbanc@in.tum.de>
parents: 784
diff changeset
   467
             val rtrm' = #rconst (qconsts_lookup thy qtrm) handle NotFound => raise exc1
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   468
           in 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   469
             if Pattern.matches thy (rtrm', rtrm) 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   470
             then rtrm else raise exc2
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   471
           end
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   472
       end 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   473
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   474
  | (t1 $ t2, t1' $ t2') =>
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   475
       (regularize_trm ctxt (t1, t1')) $ (regularize_trm ctxt (t2, t2'))
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   476
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   477
  | (Bound i, Bound i') =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   478
       if i = i' then rtrm 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   479
       else raise (LIFT_MATCH "regularize (bounds mismatch)")
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   480
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   481
  | _ =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   482
       let 
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   483
         val rtrm_str = Syntax.string_of_term ctxt rtrm
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   484
         val qtrm_str = Syntax.string_of_term ctxt qtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   485
       in
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   486
         raise (LIFT_MATCH ("regularize failed (default: " ^ rtrm_str ^ "," ^ qtrm_str ^ ")"))
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   487
       end
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   488
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   489
fun regularize_trm_chk ctxt (rtrm, qtrm) =
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   490
  regularize_trm ctxt (rtrm, qtrm) 
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   491
  |> Syntax.check_term ctxt
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   492
797
35436401f00d added a functor that allows checking what is added to the theorem lists
Christian Urban <urbanc@in.tum.de>
parents: 796
diff changeset
   493
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   494
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   495
(*** Rep/Abs Injection ***)
795
a28f805df355 renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy
Christian Urban <urbanc@in.tum.de>
parents: 792
diff changeset
   496
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   497
(*
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   498
Injection of Rep/Abs means:
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   499
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   500
  For abstractions:
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   501
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   502
  * If the type of the abstraction needs lifting, then we add Rep/Abs 
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   503
    around the abstraction; otherwise we leave it unchanged.
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   504
 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   505
  For applications:
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   506
  
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   507
  * If the application involves a bounded quantifier, we recurse on 
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   508
    the second argument. If the application is a bounded abstraction,
782
86c7ed9f354f cleaed a bit function mk_typedef_main
Christian Urban <urbanc@in.tum.de>
parents: 779
diff changeset
   509
    we always put an Rep/Abs around it (since bounded abstractions
86c7ed9f354f cleaed a bit function mk_typedef_main
Christian Urban <urbanc@in.tum.de>
parents: 779
diff changeset
   510
    are assumed to always need lifting). Otherwise we recurse on both 
86c7ed9f354f cleaed a bit function mk_typedef_main
Christian Urban <urbanc@in.tum.de>
parents: 779
diff changeset
   511
    arguments.
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   512
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   513
  For constants:
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   514
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   515
  * If the constant is (op =), we leave it always unchanged. 
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   516
    Otherwise the type of the constant needs lifting, we put
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   517
    and Rep/Abs around it. 
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   518
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   519
  For free variables:
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   520
797
35436401f00d added a functor that allows checking what is added to the theorem lists
Christian Urban <urbanc@in.tum.de>
parents: 796
diff changeset
   521
  * We put a Rep/Abs around it if the type needs lifting.
760
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   522
c1989de100b4 various tunings; map_lookup now raises an exception; addition to FIXME-TODO
Christian Urban <urbanc@in.tum.de>
parents: 758
diff changeset
   523
  Vars case cannot occur.
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   524
*)
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   525
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   526
fun mk_repabs ctxt (T, T') trm = 
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   527
  absrep_fun repF ctxt (T, T') $ (absrep_fun absF ctxt (T, T') $ trm)
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   528
833
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   529
fun inj_repabs_err ctxt msg rtrm qtrm =
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   530
let
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   531
  val rtrm_str = Syntax.string_of_term ctxt rtrm
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   532
  val qtrm_str = Syntax.string_of_term ctxt qtrm 
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   533
in
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   534
  raise LIFT_MATCH (space_implode " " [msg, quote rtrm_str, "and", quote qtrm_str])
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   535
end
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   536
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   537
849
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   538
(* bound variables need to be treated properly,
fa2b4b7af755 modifying comments/indentation in quotient_term.ml
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents: 836
diff changeset
   539
   as the type of subterms needs to be calculated   *)
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   540
fun inj_repabs_trm ctxt (rtrm, qtrm) =
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   541
 case (rtrm, qtrm) of
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   542
    (Const (@{const_name "Ball"}, T) $ r $ t, Const (@{const_name "All"}, _) $ t') =>
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   543
       Const (@{const_name "Ball"}, T) $ r $ (inj_repabs_trm ctxt (t, t'))
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   544
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   545
  | (Const (@{const_name "Bex"}, T) $ r $ t, Const (@{const_name "Ex"}, _) $ t') =>
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   546
       Const (@{const_name "Bex"}, T) $ r $ (inj_repabs_trm ctxt (t, t'))
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   547
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   548
  | (Const (@{const_name "Babs"}, T) $ r $ t, t' as (Abs _)) =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   549
      let
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   550
        val rty = fastype_of rtrm
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   551
        val qty = fastype_of qtrm
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   552
      in
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   553
        mk_repabs ctxt (rty, qty) (Const (@{const_name "Babs"}, T) $ r $ (inj_repabs_trm ctxt (t, t')))
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   554
      end
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   555
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   556
  | (Abs (x, T, t), Abs (x', T', t')) =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   557
      let
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   558
        val rty = fastype_of rtrm
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   559
        val qty = fastype_of qtrm
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   560
        val (y, s) = Term.dest_abs (x, T, t)
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   561
        val (_, s') = Term.dest_abs (x', T', t')
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   562
        val yvar = Free (y, T)
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   563
        val result = Term.lambda_name (y, yvar) (inj_repabs_trm ctxt (s, s'))
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   564
      in
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   565
        if rty = qty then result
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   566
        else mk_repabs ctxt (rty, qty) result
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   567
      end
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   568
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   569
  | (t $ s, t' $ s') =>  
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   570
       (inj_repabs_trm ctxt (t, t')) $ (inj_repabs_trm ctxt (s, s'))
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   571
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   572
  | (Free (_, T), Free (_, T')) => 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   573
        if T = T' then rtrm 
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   574
        else mk_repabs ctxt (T, T') rtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   575
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   576
  | (_, Const (@{const_name "op ="}, _)) => rtrm
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   577
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   578
  | (_, Const (_, T')) =>
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   579
      let
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   580
        val rty = fastype_of rtrm
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   581
      in 
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   582
        if rty = T' then rtrm
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   583
        else mk_repabs ctxt (rty, T') rtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   584
      end   
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   585
  
833
129caba33c03 the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
Christian Urban <urbanc@in.tum.de>
parents: 832
diff changeset
   586
  | _ => inj_repabs_err ctxt "injection (default):" rtrm qtrm
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   587
779
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   588
fun inj_repabs_trm_chk ctxt (rtrm, qtrm) =
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   589
  inj_repabs_trm ctxt (rtrm, qtrm) 
3b21b24a5fb6 corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file
Christian Urban <urbanc@in.tum.de>
parents: 776
diff changeset
   590
  |> Syntax.check_term ctxt
776
d1064fa29424 renamed get_fun to absrep_fun; introduced explicit checked versions of the term functions
Christian Urban <urbanc@in.tum.de>
parents: 775
diff changeset
   591
758
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   592
end; (* structure *)
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   593
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   594
3104d62e7a16 moved the QuotMain code into two ML-files
Christian Urban <urbanc@in.tum.de>
parents:
diff changeset
   595