| author | wenzelm | 
| Fri, 09 Jul 2021 14:41:22 +0200 | |
| changeset 73953 | 0b5e6851c722 | 
| parent 73031 | f93f0597f4fb | 
| child 74121 | bc03b0b82fe6 | 
| permissions | -rw-r--r-- | 
| 43730 | 1 | /* Title: Pure/term.scala | 
| 2 | Author: Makarius | |
| 3 | ||
| 43779 | 4 | Lambda terms, types, sorts. | 
| 43730 | 5 | |
| 6 | Note: Isabelle/ML is the primary environment for logical operations. | |
| 7 | */ | |
| 8 | ||
| 9 | package isabelle | |
| 10 | ||
| 11 | ||
| 12 | object Term | |
| 13 | {
 | |
| 70383 
38ac2e714729
more operations (avoid clones in Isabelle/MMT and Isabelle/Dedukti);
 wenzelm parents: 
68265diff
changeset | 14 | /* types and terms */ | 
| 
38ac2e714729
more operations (avoid clones in Isabelle/MMT and Isabelle/Dedukti);
 wenzelm parents: 
68265diff
changeset | 15 | |
| 70852 | 16 | sealed case class Indexname(name: String, index: Int = 0) | 
| 70537 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 17 |   {
 | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 18 | override def toString: String = | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 19 | if (index == -1) name | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 20 |       else {
 | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 21 | val dot = | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 22 |           Symbol.explode(name).reverse match {
 | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 23 | case _ :: s :: _ if s == Symbol.sub_decoded || s == Symbol.sub => false | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 24 | case c :: _ => Symbol.is_digit(c) | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 25 | case _ => true | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 26 | } | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 27 | if (dot) "?" + name + "." + index | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 28 | else if (index != 0) "?" + name + index | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 29 | else "?" + name | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 30 | } | 
| 
17160e0a60b6
Indexname.toString according to string_of_vname' in ML;
 wenzelm parents: 
70536diff
changeset | 31 | } | 
| 43730 | 32 | |
| 70850 | 33 | type Class = String | 
| 34 | type Sort = List[Class] | |
| 43730 | 35 | |
| 36 | sealed abstract class Typ | |
| 37 | case class Type(name: String, args: List[Typ] = Nil) extends Typ | |
| 70846 | 38 |   {
 | 
| 39 | override def toString: String = | |
| 40 | if (this == dummyT) "_" | |
| 41 |       else "Type(" + name + (if (args.isEmpty) "" else "," + args) + ")"
 | |
| 42 | } | |
| 70851 | 43 | case class TFree(name: String, sort: Sort = Nil) extends Typ | 
| 70846 | 44 |   {
 | 
| 45 | override def toString: String = | |
| 70851 | 46 |       "TFree(" + name + (if (sort.isEmpty) "" else "," + sort) + ")"
 | 
| 70846 | 47 | } | 
| 70851 | 48 | case class TVar(name: Indexname, sort: Sort = Nil) extends Typ | 
| 70846 | 49 |   {
 | 
| 50 | override def toString: String = | |
| 70851 | 51 |       "TVar(" + name + (if (sort.isEmpty) "" else "," + sort) + ")"
 | 
| 70846 | 52 | } | 
| 71601 | 53 |   val dummyT: Type = Type("dummy")
 | 
| 43730 | 54 | |
| 55 | sealed abstract class Term | |
| 71221 | 56 |   {
 | 
| 57 | def head: Term = | |
| 58 |       this match {
 | |
| 59 | case App(fun, _) => fun.head | |
| 60 | case _ => this | |
| 61 | } | |
| 62 | } | |
| 70846 | 63 | case class Const(name: String, typargs: List[Typ] = Nil) extends Term | 
| 64 |   {
 | |
| 65 | override def toString: String = | |
| 70897 | 66 | if (this == dummy) "_" | 
| 67 |       else "Const(" + name + (if (typargs.isEmpty) "" else "," + typargs) + ")"
 | |
| 70846 | 68 | } | 
| 43730 | 69 | case class Free(name: String, typ: Typ = dummyT) extends Term | 
| 70846 | 70 |   {
 | 
| 71 | override def toString: String = | |
| 72 |       "Free(" + name + (if (typ == dummyT) "" else "," + typ) + ")"
 | |
| 73 | } | |
| 43730 | 74 | case class Var(name: Indexname, typ: Typ = dummyT) extends Term | 
| 70846 | 75 |   {
 | 
| 76 | override def toString: String = | |
| 77 |       "Var(" + name + (if (typ == dummyT) "" else "," + typ) + ")"
 | |
| 78 | } | |
| 43730 | 79 | case class Bound(index: Int) extends Term | 
| 70846 | 80 | case class Abs(name: String, typ: Typ, body: Term) extends Term | 
| 43730 | 81 | case class App(fun: Term, arg: Term) extends Term | 
| 70850 | 82 |   {
 | 
| 83 | override def toString: String = | |
| 84 |       this match {
 | |
| 85 |         case OFCLASS(ty, c) => "OFCLASS(" + ty + "," + c + ")"
 | |
| 86 |         case _ => "App(" + fun + "," + arg + ")"
 | |
| 87 | } | |
| 88 | } | |
| 68265 | 89 | |
| 70897 | 90 |   def dummy_pattern(ty: Typ): Term = Const("Pure.dummy_pattern", List(ty))
 | 
| 91 | val dummy: Term = dummy_pattern(dummyT) | |
| 92 | ||
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 93 | sealed abstract class Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 94 | case object MinProof extends Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 95 | case class PBound(index: Int) extends Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 96 | case class Abst(name: String, typ: Typ, body: Proof) extends Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 97 | case class AbsP(name: String, hyp: Term, body: Proof) extends Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 98 | case class Appt(fun: Proof, arg: Term) extends Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 99 | case class AppP(fun: Proof, arg: Proof) extends Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 100 | case class Hyp(hyp: Term) extends Proof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 101 | case class PAxm(name: String, types: List[Typ]) extends Proof | 
| 71777 
3875815f5967
clarified signature: avoid clash with Isabelle/Scala Term.OFCLASS on case-insensible file-system;
 wenzelm parents: 
71601diff
changeset | 102 | case class PClass(typ: Typ, cls: Class) extends Proof | 
| 70834 | 103 | case class Oracle(name: String, prop: Term, types: List[Typ]) extends Proof | 
| 70916 
4c15217d6266
clarified signature: name of standard_proof is authentic, otherwise empty;
 wenzelm parents: 
70897diff
changeset | 104 | case class PThm(serial: Long, theory_name: String, name: String, types: List[Typ]) extends Proof | 
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 105 | |
| 68265 | 106 | |
| 70850 | 107 | /* type classes within the logic */ | 
| 70385 
68d2c533db9c
more operations: support type classes within the logic;
 wenzelm parents: 
70383diff
changeset | 108 | |
| 70850 | 109 | object Class_Const | 
| 110 |   {
 | |
| 111 | val suffix = "_class" | |
| 112 | def apply(c: Class): String = c + suffix | |
| 113 | def unapply(s: String): Option[Class] = | |
| 114 | if (s.endsWith(suffix)) Some(s.substring(0, s.length - suffix.length)) else None | |
| 115 | } | |
| 70385 
68d2c533db9c
more operations: support type classes within the logic;
 wenzelm parents: 
70383diff
changeset | 116 | |
| 70850 | 117 | object OFCLASS | 
| 118 |   {
 | |
| 119 | def apply(ty: Typ, s: Sort): List[Term] = s.map(c => apply(ty, c)) | |
| 120 | ||
| 121 | def apply(ty: Typ, c: Class): Term = | |
| 122 | App(Const(Class_Const(c), List(ty)), Const(Pure_Thy.TYPE, List(ty))) | |
| 70385 
68d2c533db9c
more operations: support type classes within the logic;
 wenzelm parents: 
70383diff
changeset | 123 | |
| 70850 | 124 | def unapply(t: Term): Option[(Typ, String)] = | 
| 125 |       t match {
 | |
| 126 | case App(Const(Class_Const(c), List(ty)), Const(Pure_Thy.TYPE, List(ty1))) | |
| 127 | if ty == ty1 => Some((ty, c)) | |
| 128 | case _ => None | |
| 129 | } | |
| 70385 
68d2c533db9c
more operations: support type classes within the logic;
 wenzelm parents: 
70383diff
changeset | 130 | } | 
| 
68d2c533db9c
more operations: support type classes within the logic;
 wenzelm parents: 
70383diff
changeset | 131 | |
| 
68d2c533db9c
more operations: support type classes within the logic;
 wenzelm parents: 
70383diff
changeset | 132 | |
| 68265 | 133 | |
| 134 | /** cache **/ | |
| 135 | ||
| 73024 | 136 | object Cache | 
| 137 |   {
 | |
| 138 | def make( | |
| 73026 
237bd6318cc1
more uniform default --- hardly relevant in practice;
 wenzelm parents: 
73024diff
changeset | 139 | max_string: Int = isabelle.Cache.default_max_string, | 
| 73024 | 140 | initial_size: Int = isabelle.Cache.default_initial_size): Cache = | 
| 141 | new Cache(initial_size, max_string) | |
| 68265 | 142 | |
| 73024 | 143 | val none: Cache = make(max_string = 0) | 
| 144 | } | |
| 145 | ||
| 146 | class Cache private[Term](max_string: Int, initial_size: Int) | |
| 73031 
f93f0597f4fb
clarified signature: absorb XZ.Cache into XML.Cache;
 wenzelm parents: 
73026diff
changeset | 147 | extends isabelle.Cache(max_string, initial_size) | 
| 68265 | 148 |   {
 | 
| 149 | protected def cache_indexname(x: Indexname): Indexname = | |
| 70536 | 150 | lookup(x) getOrElse store(Indexname(cache_string(x.name), x.index)) | 
| 68265 | 151 | |
| 152 | protected def cache_sort(x: Sort): Sort = | |
| 73024 | 153 | if (x.isEmpty) Nil | 
| 154 | else lookup(x) getOrElse store(x.map(cache_string)) | |
| 68265 | 155 | |
| 156 | protected def cache_typ(x: Typ): Typ = | |
| 157 |     {
 | |
| 158 | if (x == dummyT) dummyT | |
| 159 | else | |
| 160 |         lookup(x) match {
 | |
| 161 | case Some(y) => y | |
| 162 | case None => | |
| 163 |             x match {
 | |
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 164 | case Type(name, args) => store(Type(cache_string(name), cache_typs(args))) | 
| 68265 | 165 | case TFree(name, sort) => store(TFree(cache_string(name), cache_sort(sort))) | 
| 166 | case TVar(name, sort) => store(TVar(cache_indexname(name), cache_sort(sort))) | |
| 167 | } | |
| 168 | } | |
| 169 | } | |
| 170 | ||
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 171 | protected def cache_typs(x: List[Typ]): List[Typ] = | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 172 |     {
 | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 173 | if (x.isEmpty) Nil | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 174 |       else {
 | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 175 |         lookup(x) match {
 | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 176 | case Some(y) => y | 
| 71601 | 177 | case None => store(x.map(cache_typ)) | 
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 178 | } | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 179 | } | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 180 | } | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 181 | |
| 68265 | 182 | protected def cache_term(x: Term): Term = | 
| 183 |     {
 | |
| 184 |       lookup(x) match {
 | |
| 185 | case Some(y) => y | |
| 186 | case None => | |
| 187 |           x match {
 | |
| 70784 
799437173553
Term_XML.Encode/Decode.term uses Const "typargs";
 wenzelm parents: 
70559diff
changeset | 188 | case Const(name, typargs) => store(Const(cache_string(name), cache_typs(typargs))) | 
| 68265 | 189 | case Free(name, typ) => store(Free(cache_string(name), cache_typ(typ))) | 
| 190 | case Var(name, typ) => store(Var(cache_indexname(name), cache_typ(typ))) | |
| 70536 | 191 | case Bound(_) => store(x) | 
| 68265 | 192 | case Abs(name, typ, body) => | 
| 193 | store(Abs(cache_string(name), cache_typ(typ), cache_term(body))) | |
| 194 | case App(fun, arg) => store(App(cache_term(fun), cache_term(arg))) | |
| 195 | } | |
| 196 | } | |
| 197 | } | |
| 198 | ||
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 199 | protected def cache_proof(x: Proof): Proof = | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 200 |     {
 | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 201 | if (x == MinProof) MinProof | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 202 |       else {
 | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 203 |         lookup(x) match {
 | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 204 | case Some(y) => y | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 205 | case None => | 
| 71781 | 206 |             (x: @unchecked) match {
 | 
| 70536 | 207 | case PBound(_) => store(x) | 
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 208 | case Abst(name, typ, body) => | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 209 | store(Abst(cache_string(name), cache_typ(typ), cache_proof(body))) | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 210 | case AbsP(name, hyp, body) => | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 211 | store(AbsP(cache_string(name), cache_term(hyp), cache_proof(body))) | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 212 | case Appt(fun, arg) => store(Appt(cache_proof(fun), cache_term(arg))) | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 213 | case AppP(fun, arg) => store(AppP(cache_proof(fun), cache_proof(arg))) | 
| 70535 | 214 | case Hyp(hyp) => store(Hyp(cache_term(hyp))) | 
| 215 | case PAxm(name, types) => store(PAxm(cache_string(name), cache_typs(types))) | |
| 71777 
3875815f5967
clarified signature: avoid clash with Isabelle/Scala Term.OFCLASS on case-insensible file-system;
 wenzelm parents: 
71601diff
changeset | 216 | case PClass(typ, cls) => store(PClass(cache_typ(typ), cache_string(cls))) | 
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 217 | case Oracle(name, prop, types) => | 
| 70834 | 218 | store(Oracle(cache_string(name), cache_term(prop), cache_typs(types))) | 
| 70538 
fc9ba6fe367f
clarified PThm: theory_name simplifies retrieval from exports;
 wenzelm parents: 
70537diff
changeset | 219 | case PThm(serial, theory_name, name, types) => | 
| 
fc9ba6fe367f
clarified PThm: theory_name simplifies retrieval from exports;
 wenzelm parents: 
70537diff
changeset | 220 | store(PThm(serial, cache_string(theory_name), cache_string(name), cache_typs(types))) | 
| 70533 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 221 | } | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 222 | } | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 223 | } | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 224 | } | 
| 
031620901fcd
support for (fully reconstructed) proof terms in Scala;
 wenzelm parents: 
70385diff
changeset | 225 | |
| 68265 | 226 | // main methods | 
| 73024 | 227 | def indexname(x: Indexname): Indexname = | 
| 228 |       if (no_cache) x else synchronized { cache_indexname(x) }
 | |
| 229 | def sort(x: Sort): Sort = | |
| 230 |       if (no_cache) x else synchronized { cache_sort(x) }
 | |
| 231 | def typ(x: Typ): Typ = | |
| 232 |       if (no_cache) x else synchronized { cache_typ(x) }
 | |
| 233 | def term(x: Term): Term = | |
| 234 |       if (no_cache) x else synchronized { cache_term(x) }
 | |
| 235 | def proof(x: Proof): Proof = | |
| 236 |       if (no_cache) x else synchronized { cache_proof(x) }
 | |
| 68265 | 237 | |
| 238 | def position(x: Position.T): Position.T = | |
| 73024 | 239 | if (no_cache) x | 
| 240 |       else synchronized { x.map({ case (a, b) => (cache_string(a), cache_string(b)) }) }
 | |
| 68265 | 241 | } | 
| 43731 
70072780e095
inner syntax supports inlined YXML according to Term_XML (particularly useful for producing text under program control);
 wenzelm parents: 
43730diff
changeset | 242 | } |